Skip to content

Commit

Permalink
Only export R from Rbase to avoid name clashes
Browse files Browse the repository at this point in the history
In particular, there's a constructor called IRQ.
  • Loading branch information
bacam committed Nov 14, 2023
1 parent c20045e commit fa0c524
Showing 1 changed file with 3 additions and 1 deletion.
4 changes: 3 additions & 1 deletion src/Real.v
Original file line number Diff line number Diff line change
Expand Up @@ -65,13 +65,15 @@
(* SUCH DAMAGE. *)
(*==========================================================================*)

Require Export Rbase.
Require Import Rbase.
Require Import Reals.
Require Export ROrderedType.
Require Import Sail.Values.
Require Import Lia.
Local Open Scope Z.

Export Rdefinitions(R).

(* "Decidable" in a classical sense... *)
#[export] Instance Decidable_eq_real : forall (x y : R), Decidable (x = y) :=
Decidable_eq_from_dec Req_dec.
Expand Down

0 comments on commit fa0c524

Please sign in to comment.