Skip to content
Open
Show file tree
Hide file tree
Changes from all commits
Commits
File filter

Filter by extension

Filter by extension

Conversations
Failed to load comments.
Loading
Jump to
Jump to file
Failed to load files.
Loading
Diff view
Diff view
4 changes: 2 additions & 2 deletions theories/cauchyreals.v
Original file line number Diff line number Diff line change
Expand Up @@ -628,7 +628,7 @@ Lemma cst_crealP (x : F) : creal_axiom (fun _ => x).
Proof. by exists (fun _ => 0%N)=> *; rewrite subrr normr0. Qed.
Definition cst_creal (x : F) := CReal (cst_crealP x).
Notation "x %:CR" := (cst_creal x)
(at level 2, left associativity, format "x %:CR") : creal_scope.
(at level 1, left associativity, format "x %:CR") : creal_scope.
Notation "0" := (0 %:CR) : creal_scope.

Lemma lbound0P (x : creal) (x_neq0 : x != 0) i :
Expand Down Expand Up @@ -1638,7 +1638,7 @@ Notation "!=%CR" := neq_creal : creal_scope.
Notation "x != y" := (neq_creal x y) : creal_scope.

Notation "x %:CR" := (cst_creal x)
(at level 2, left associativity, format "x %:CR") : creal_scope.
(at level 1, left associativity, format "x %:CR") : creal_scope.
Notation "0" := (0 %:CR)%CR : creal_scope.

Notation "<%CR" := lt_creal : creal_scope.
Expand Down
2 changes: 1 addition & 1 deletion theories/complex.v
Original file line number Diff line number Diff line change
Expand Up @@ -30,7 +30,7 @@ Reserved Notation "x +i* y"
Reserved Notation "x -i* y"
(at level 40, left associativity, format "x -i* y").
Reserved Notation "R [i]"
(at level 2, left associativity, format "R [i]").
(at level 1, left associativity, format "R [i]").

Local Notation sgr := Num.sg.
Local Notation sqrtr := Num.sqrt.
Expand Down
6 changes: 3 additions & 3 deletions theories/realalg.v
Original file line number Diff line number Diff line change
Expand Up @@ -571,7 +571,7 @@ Definition to_alg_def (phF : phant F) : F -> alg :=
lift_embed alg cst_algcreal.
Notation to_alg := (@to_alg_def (Phant F)).
Notation "x %:RA" := (to_alg x)
(at level 2, left associativity, format "x %:RA").
(at level 1, left associativity, format "x %:RA").
Local Notation "p ^ f" := (map_poly f p) : ring_scope.

Canonical to_alg_pi_morph := PiEmbed to_alg.
Expand Down Expand Up @@ -1176,7 +1176,7 @@ End RealAlg.

Notation to_alg F := (@to_alg_def _ (Phant F)).
Notation "x %:RA" := (to_alg _ x)
(at level 2, left associativity, format "x %:RA").
(at level 1, left associativity, format "x %:RA").

Lemma upper_nthrootVP (F : archiFieldType) (x : F) (i : nat) :
0 < x -> (Num.bound (x ^-1) <= i)%N -> 2%:R ^- i < x.
Expand Down Expand Up @@ -1381,7 +1381,7 @@ Notation "{ 'realclosure' F }" := (RealAlg.alg F).
Notation annul_realalg := RealAlg.annul_alg.
Notation realalg_of F := (@RealAlg.to_alg_def _ (Phant F)).
Notation "x %:RA" := (realalg_of x)
(at level 2, left associativity, format "x %:RA").
(at level 1, left associativity, format "x %:RA").

HB.instance Definition _ (F : archiFieldType) := GRing.RMorphism.on (to_alg F).

Expand Down