We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent f39bbcf commit 5435910Copy full SHA for 5435910
Cslib/Foundations/Semantics/LTS/Bisimulation.lean
@@ -235,11 +235,11 @@ section Order
235
236
/-! ## Order properties -/
237
238
-noncomputable instance : Max {r // lts.IsBisimulation r} where
+instance : Max {r // lts.IsBisimulation r} where
239
max r s := ⟨r.1 ⊔ s.1, Bisimulation.union r.2 s.2⟩
240
241
/-- Bisimulations equipped with union form a join-semilattice. -/
242
-noncomputable instance : SemilatticeSup {r // lts.IsBisimulation r} where
+instance : SemilatticeSup {r // lts.IsBisimulation r} where
243
sup r s := r ⊔ s
244
le_sup_left r s := by
245
simp only [LE.le]
0 commit comments