Skip to content

Commit

Permalink
Merge pull request #129 from leanprover-community/more_example_updates
Browse files Browse the repository at this point in the history
  • Loading branch information
jcommelin committed Oct 14, 2022
2 parents ebb498c + bdb33ea commit 92f188b
Show file tree
Hide file tree
Showing 3 changed files with 5 additions and 5 deletions.
2 changes: 1 addition & 1 deletion src/examples/Ext.lean
Expand Up @@ -92,7 +92,7 @@ rfl
`Ext' 0 (X, Y) β‰… Hom(X,Y)`.
-/
example (X Y : 𝓐) : Ext' 0 (op X) Y β‰… AddCommGroup.of (X ⟢ Y) :=
(Ext'_zero_flip_iso _ _).app _
(Ext'_zero_flip_iso 𝓐 Y).app (op X)

/-!
The isomorphism above is functorial in the first variable, and the isomorphism of functors
Expand Down
4 changes: 2 additions & 2 deletions src/examples/cond.lean
Expand Up @@ -118,8 +118,8 @@ example
(Ο€ : Ξ  i, X i ⟢ B)
-- such that `Ο€` is jointly surjective,
(hΟ€ : βˆ€ b : B, βˆƒ i (x : X i), Ο€ i x = b)
-- and all families of elements `x i : F (op $ X i)`,
(x : Ξ  i, F (op $ X i))
-- and all families of elements `x i : F (op (X i))`,
(x : Ξ  i, F (op (X i)))
-- which are compatible on pullbacks `X i Γ—_{B} X j`
(hx : βˆ€ i j : Ξ±,
F.map (pullback.fst : pullback (Ο€ i) (Ο€ j) ⟢ X i).op (x i) =
Expand Down
4 changes: 2 additions & 2 deletions src/examples/real.lean
Expand Up @@ -32,12 +32,12 @@ rfl
/-!
Any conditionally complete linear ordered field is isomorphic (as an ordered ring) to `ℝ`.
-/
example {R : Type*} [conditionally_complete_linear_ordered_field R] : R ≃+*o ℝ :=
example {R : Type} [conditionally_complete_linear_ordered_field R] : R ≃+*o ℝ :=
default

/-!
The isomorphism above is unique.
-/
example {R : Type*} [conditionally_complete_linear_ordered_field R] (e₁ eβ‚‚ : R ≃+*o ℝ) :
example {R : Type} [conditionally_complete_linear_ordered_field R] (e₁ eβ‚‚ : R ≃+*o ℝ) :
e₁ = eβ‚‚ :=
subsingleton.elim _ _

0 comments on commit 92f188b

Please sign in to comment.