src/HOLCF/domain/axioms.ML
author wenzelm
Thu, 14 Jul 2005 19:28:24 +0200
changeset 16842 5979c46853d1
parent 16778 2162c0de4673
child 17811 10ebcd7032c1
permissions -rw-r--r--
tuned;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
2453
2d416226b27d corrected headers
oheimb
parents: 1637
diff changeset
     1
(*  Title:      HOLCF/domain/axioms.ML
2d416226b27d corrected headers
oheimb
parents: 1637
diff changeset
     2
    ID:         $Id$
12030
wenzelm
parents: 11531
diff changeset
     3
    Author:     David von Oheimb
2453
2d416226b27d corrected headers
oheimb
parents: 1637
diff changeset
     4
12030
wenzelm
parents: 11531
diff changeset
     5
Syntax generator for domain section.
1274
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
     6
*)
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
     7
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
     8
structure Domain_Axioms = struct
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
     9
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    10
local
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    11
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    12
open Domain_Library;
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    13
infixr 0 ===>;infixr 0 ==>;infix 0 == ; 
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    14
infix 1 ===; infix 1 ~= ; infix 1 <<; infix 1 ~<<;
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    15
infix 9 `   ; infix 9 `% ; infix 9 `%%; infixr 9 oo;
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    16
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    17
fun infer_types thy' = map (inferT_axm (sign_of thy'));
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    18
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    19
fun calc_axioms comp_dname (eqs : eq list) n (((dname,_),cons) : eq)=
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    20
let
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    21
1637
b8a8ae2e5de1 Updated: 01-Mar-96 when functional strictified, copy_def based on when_def
oheimb
parents: 1461
diff changeset
    22
(* ----- axioms and definitions concerning the isomorphism ------------------ *)
1274
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    23
11531
d038246a62f2 Renamed functions % and %% to avoid clash with syntax for proof terms.
berghofe
parents: 8438
diff changeset
    24
  val dc_abs = %%:(dname^"_abs");
d038246a62f2 Renamed functions % and %% to avoid clash with syntax for proof terms.
berghofe
parents: 8438
diff changeset
    25
  val dc_rep = %%:(dname^"_rep");
1274
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    26
  val x_name'= "x";
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    27
  val x_name = idx_name eqs x_name' (n+1);
4008
2444085532c6 adapted domain and ax_ops package for name spaces
oheimb
parents: 3771
diff changeset
    28
  val dnam = Sign.base_name dname;
1274
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    29
11531
d038246a62f2 Renamed functions % and %% to avoid clash with syntax for proof terms.
berghofe
parents: 8438
diff changeset
    30
 val abs_iso_ax = ("abs_iso" ,mk_trp(dc_rep`(dc_abs`%x_name')=== %:x_name'));
d038246a62f2 Renamed functions % and %% to avoid clash with syntax for proof terms.
berghofe
parents: 8438
diff changeset
    31
 val rep_iso_ax = ("rep_iso" ,mk_trp(dc_abs`(dc_rep`%x_name')=== %:x_name'));
1274
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    32
11531
d038246a62f2 Renamed functions % and %% to avoid clash with syntax for proof terms.
berghofe
parents: 8438
diff changeset
    33
  val when_def = ("when_def",%%:(dname^"_when") == 
15574
b1d1b5bfc464 Removed practically all references to Library.foldr.
skalberg
parents: 15570
diff changeset
    34
     foldr (uncurry /\ ) (/\x_name'((when_body cons (fn (x,y) =>
b1d1b5bfc464 Removed practically all references to Library.foldr.
skalberg
parents: 15570
diff changeset
    35
				Bound(1+length cons+x-y)))`(dc_rep`Bound 0))) (when_funs cons));
1274
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    36
1637
b8a8ae2e5de1 Updated: 01-Mar-96 when functional strictified, copy_def based on when_def
oheimb
parents: 1461
diff changeset
    37
  fun con_def outer recu m n (_,args) = let
16842
wenzelm
parents: 16778
diff changeset
    38
     fun idxs z x arg = (if is_lazy arg then fn t => %%:upN`t else I)
4755
843b5f159c7e added cproj', and therefore extended prj
oheimb
parents: 4122
diff changeset
    39
			(if recu andalso is_rec arg then (cproj (Bound z) eqs
843b5f159c7e added cproj', and therefore extended prj
oheimb
parents: 4122
diff changeset
    40
				  (rec_of arg))`Bound(z-x) else Bound(z-x));
16778
2162c0de4673 use qualified names for all constants
huffman
parents: 16394
diff changeset
    41
     fun parms [] = %%:ONE_N
2162c0de4673 use qualified names for all constants
huffman
parents: 16394
diff changeset
    42
     |   parms vs = foldr'(fn(x,t)=> %%:spairN`x`t)(mapn (idxs(length vs))1 vs);
1637
b8a8ae2e5de1 Updated: 01-Mar-96 when functional strictified, copy_def based on when_def
oheimb
parents: 1461
diff changeset
    43
     fun inj y 1 _ = y
16778
2162c0de4673 use qualified names for all constants
huffman
parents: 16394
diff changeset
    44
     |   inj y _ 0 = %%:sinlN`y
2162c0de4673 use qualified names for all constants
huffman
parents: 16394
diff changeset
    45
     |   inj y i j = %%:sinrN`(inj y (i-1) (j-1));
15574
b1d1b5bfc464 Removed practically all references to Library.foldr.
skalberg
parents: 15570
diff changeset
    46
  in foldr /\# (outer (inj (parms args) m n)) args end;
1274
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    47
11531
d038246a62f2 Renamed functions % and %% to avoid clash with syntax for proof terms.
berghofe
parents: 8438
diff changeset
    48
  val copy_def = ("copy_def", %%:(dname^"_copy") == /\"f" (dc_abs oo 
15570
8d8c70b41bab Move towards standard functions.
skalberg
parents: 14981
diff changeset
    49
	Library.foldl (op `) (%%:(dname^"_when") , 
16842
wenzelm
parents: 16778
diff changeset
    50
	              mapn (con_def I true (length cons)) 0 cons)));
1274
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    51
1637
b8a8ae2e5de1 Updated: 01-Mar-96 when functional strictified, copy_def based on when_def
oheimb
parents: 1461
diff changeset
    52
(* -- definitions concerning the constructors, discriminators and selectors - *)
b8a8ae2e5de1 Updated: 01-Mar-96 when functional strictified, copy_def based on when_def
oheimb
parents: 1461
diff changeset
    53
4043
35766855f344 domain package:
oheimb
parents: 4008
diff changeset
    54
  val con_defs = mapn (fn n => fn (con,args) => (extern_name con ^"_def",  
11531
d038246a62f2 Renamed functions % and %% to avoid clash with syntax for proof terms.
berghofe
parents: 8438
diff changeset
    55
  %%:con == con_def (fn t => dc_abs`t) false (length cons) n (con,args))) 0 cons;
1274
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    56
4043
35766855f344 domain package:
oheimb
parents: 4008
diff changeset
    57
  val dis_defs = let
11531
d038246a62f2 Renamed functions % and %% to avoid clash with syntax for proof terms.
berghofe
parents: 8438
diff changeset
    58
	fun ddef (con,_) = (dis_name con ^"_def",%%:(dis_name con) == 
d038246a62f2 Renamed functions % and %% to avoid clash with syntax for proof terms.
berghofe
parents: 8438
diff changeset
    59
		 mk_cRep_CFun(%%:(dname^"_when"),map 
15574
b1d1b5bfc464 Removed practically all references to Library.foldr.
skalberg
parents: 15570
diff changeset
    60
			(fn (con',args) => (foldr /\#
16778
2162c0de4673 use qualified names for all constants
huffman
parents: 16394
diff changeset
    61
			   (if con'=con then %%:TT_N else %%:FF_N) args)) cons))
1637
b8a8ae2e5de1 Updated: 01-Mar-96 when functional strictified, copy_def based on when_def
oheimb
parents: 1461
diff changeset
    62
	in map ddef cons end;
1274
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    63
16224
57094b83774e Domain package generates match functions for new datatypes, for use with the fixrec package
huffman
parents: 15574
diff changeset
    64
  val mat_defs = let
57094b83774e Domain package generates match functions for new datatypes, for use with the fixrec package
huffman
parents: 15574
diff changeset
    65
	fun mdef (con,_) = (mat_name con ^"_def",%%:(mat_name con) == 
57094b83774e Domain package generates match functions for new datatypes, for use with the fixrec package
huffman
parents: 15574
diff changeset
    66
		 mk_cRep_CFun(%%:(dname^"_when"),map 
57094b83774e Domain package generates match functions for new datatypes, for use with the fixrec package
huffman
parents: 15574
diff changeset
    67
			(fn (con',args) => (foldr /\#
16778
2162c0de4673 use qualified names for all constants
huffman
parents: 16394
diff changeset
    68
			   (if con'=con
2162c0de4673 use qualified names for all constants
huffman
parents: 16394
diff changeset
    69
                               then %%:returnN`(mk_ctuple (map (bound_arg args) args))
2162c0de4673 use qualified names for all constants
huffman
parents: 16394
diff changeset
    70
                               else %%:failN) args)) cons))
16224
57094b83774e Domain package generates match functions for new datatypes, for use with the fixrec package
huffman
parents: 15574
diff changeset
    71
	in map mdef cons end;
57094b83774e Domain package generates match functions for new datatypes, for use with the fixrec package
huffman
parents: 15574
diff changeset
    72
4043
35766855f344 domain package:
oheimb
parents: 4008
diff changeset
    73
  val sel_defs = let
16394
495dbcd4f4c9 in domain declarations, selector names are now optional
huffman
parents: 16332
diff changeset
    74
	fun sdef con n arg = Option.map (fn sel => (sel^"_def",%%:sel == 
11531
d038246a62f2 Renamed functions % and %% to avoid clash with syntax for proof terms.
berghofe
parents: 8438
diff changeset
    75
		 mk_cRep_CFun(%%:(dname^"_when"),map 
16778
2162c0de4673 use qualified names for all constants
huffman
parents: 16394
diff changeset
    76
			(fn (con',args) => if con'<>con then UU else
16394
495dbcd4f4c9 in domain declarations, selector names are now optional
huffman
parents: 16332
diff changeset
    77
			 foldr /\# (Bound (length args - n)) args) cons))) (sel_of arg);
16842
wenzelm
parents: 16778
diff changeset
    78
	in List.mapPartial I (List.concat(map (fn (con,args) => mapn (sdef con) 1 args) cons)) end;
1274
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    79
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    80
1637
b8a8ae2e5de1 Updated: 01-Mar-96 when functional strictified, copy_def based on when_def
oheimb
parents: 1461
diff changeset
    81
(* ----- axiom and definitions concerning induction ------------------------- *)
1274
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    82
16778
2162c0de4673 use qualified names for all constants
huffman
parents: 16394
diff changeset
    83
  val reach_ax = ("reach", mk_trp(cproj (%%:fixN`%%(comp_dname^"_copy")) eqs n
11531
d038246a62f2 Renamed functions % and %% to avoid clash with syntax for proof terms.
berghofe
parents: 8438
diff changeset
    84
					`%x_name === %:x_name));
d038246a62f2 Renamed functions % and %% to avoid clash with syntax for proof terms.
berghofe
parents: 8438
diff changeset
    85
  val take_def = ("take_def",%%:(dname^"_take") == mk_lam("n",cproj' 
16778
2162c0de4673 use qualified names for all constants
huffman
parents: 16394
diff changeset
    86
	     (%%:iterateN $ Bound 0 $ %%:(comp_dname^"_copy") $ UU) eqs n));
11531
d038246a62f2 Renamed functions % and %% to avoid clash with syntax for proof terms.
berghofe
parents: 8438
diff changeset
    87
  val finite_def = ("finite_def",%%:(dname^"_finite") == mk_lam(x_name,
d038246a62f2 Renamed functions % and %% to avoid clash with syntax for proof terms.
berghofe
parents: 8438
diff changeset
    88
	mk_ex("n",(%%:(dname^"_take") $ Bound 0)`Bound 1 === Bound 1)));
1274
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    89
4043
35766855f344 domain package:
oheimb
parents: 4008
diff changeset
    90
in (dnam,
35766855f344 domain package:
oheimb
parents: 4008
diff changeset
    91
    [abs_iso_ax, rep_iso_ax, reach_ax],
35766855f344 domain package:
oheimb
parents: 4008
diff changeset
    92
    [when_def, copy_def] @
16224
57094b83774e Domain package generates match functions for new datatypes, for use with the fixrec package
huffman
parents: 15574
diff changeset
    93
     con_defs @ dis_defs @ mat_defs @ sel_defs @
4043
35766855f344 domain package:
oheimb
parents: 4008
diff changeset
    94
    [take_def, finite_def])
1637
b8a8ae2e5de1 Updated: 01-Mar-96 when functional strictified, copy_def based on when_def
oheimb
parents: 1461
diff changeset
    95
end; (* let *)
1274
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    96
8438
b8389b4fca9c adapted to new PureThy.add_thms etc.;
wenzelm
parents: 6092
diff changeset
    97
fun add_axioms_i x = #1 o PureThy.add_axioms_i (map Thm.no_attributes x);
16332
25a440fe5f65 add_axioms_infer -- avoids use of stale theory;
wenzelm
parents: 16224
diff changeset
    98
fun add_axioms_infer axms thy = add_axioms_i (infer_types thy axms) thy;
1274
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
    99
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
   100
in (* local *)
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
   101
4008
2444085532c6 adapted domain and ax_ops package for name spaces
oheimb
parents: 3771
diff changeset
   102
fun add_axioms (comp_dnam, eqs : eq list) thy' = let
2444085532c6 adapted domain and ax_ops package for name spaces
oheimb
parents: 3771
diff changeset
   103
  val comp_dname = Sign.full_name (sign_of thy') comp_dnam;
1274
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
   104
  val dnames = map (fst o fst) eqs;
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
   105
  val x_name = idx_name dnames "x"; 
11531
d038246a62f2 Renamed functions % and %% to avoid clash with syntax for proof terms.
berghofe
parents: 8438
diff changeset
   106
  fun copy_app dname = %%:(dname^"_copy")`Bound 0;
d038246a62f2 Renamed functions % and %% to avoid clash with syntax for proof terms.
berghofe
parents: 8438
diff changeset
   107
  val copy_def = ("copy_def" , %%:(comp_dname^"_copy") ==
1637
b8a8ae2e5de1 Updated: 01-Mar-96 when functional strictified, copy_def based on when_def
oheimb
parents: 1461
diff changeset
   108
				    /\"f"(foldr' cpair (map copy_app dnames)));
11531
d038246a62f2 Renamed functions % and %% to avoid clash with syntax for proof terms.
berghofe
parents: 8438
diff changeset
   109
  val bisim_def = ("bisim_def",%%:(comp_dname^"_bisim")==mk_lam("R",
1274
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
   110
    let
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
   111
      fun one_con (con,args) = let
1637
b8a8ae2e5de1 Updated: 01-Mar-96 when functional strictified, copy_def based on when_def
oheimb
parents: 1461
diff changeset
   112
	val nonrec_args = filter_out is_rec args;
15570
8d8c70b41bab Move towards standard functions.
skalberg
parents: 14981
diff changeset
   113
	val    rec_args = List.filter     is_rec args;
1637
b8a8ae2e5de1 Updated: 01-Mar-96 when functional strictified, copy_def based on when_def
oheimb
parents: 1461
diff changeset
   114
	val    recs_cnt = length rec_args;
b8a8ae2e5de1 Updated: 01-Mar-96 when functional strictified, copy_def based on when_def
oheimb
parents: 1461
diff changeset
   115
	val allargs     = nonrec_args @ rec_args
b8a8ae2e5de1 Updated: 01-Mar-96 when functional strictified, copy_def based on when_def
oheimb
parents: 1461
diff changeset
   116
				      @ map (upd_vname (fn s=> s^"'")) rec_args;
b8a8ae2e5de1 Updated: 01-Mar-96 when functional strictified, copy_def based on when_def
oheimb
parents: 1461
diff changeset
   117
	val allvns      = map vname allargs;
b8a8ae2e5de1 Updated: 01-Mar-96 when functional strictified, copy_def based on when_def
oheimb
parents: 1461
diff changeset
   118
	fun vname_arg s arg = if is_rec arg then vname arg^s else vname arg;
b8a8ae2e5de1 Updated: 01-Mar-96 when functional strictified, copy_def based on when_def
oheimb
parents: 1461
diff changeset
   119
	val vns1        = map (vname_arg "" ) args;
b8a8ae2e5de1 Updated: 01-Mar-96 when functional strictified, copy_def based on when_def
oheimb
parents: 1461
diff changeset
   120
	val vns2        = map (vname_arg "'") args;
b8a8ae2e5de1 Updated: 01-Mar-96 when functional strictified, copy_def based on when_def
oheimb
parents: 1461
diff changeset
   121
	val allargs_cnt = length nonrec_args + 2*recs_cnt;
b8a8ae2e5de1 Updated: 01-Mar-96 when functional strictified, copy_def based on when_def
oheimb
parents: 1461
diff changeset
   122
	val rec_idxs    = (recs_cnt-1) downto 0;
b8a8ae2e5de1 Updated: 01-Mar-96 when functional strictified, copy_def based on when_def
oheimb
parents: 1461
diff changeset
   123
	val nonlazy_idxs = map snd (filter_out (fn (arg,_) => is_lazy arg)
b8a8ae2e5de1 Updated: 01-Mar-96 when functional strictified, copy_def based on when_def
oheimb
parents: 1461
diff changeset
   124
					 (allargs~~((allargs_cnt-1) downto 0)));
4755
843b5f159c7e added cproj', and therefore extended prj
oheimb
parents: 4122
diff changeset
   125
	fun rel_app i ra = proj (Bound(allargs_cnt+2)) eqs (rec_of ra) $ 
1637
b8a8ae2e5de1 Updated: 01-Mar-96 when functional strictified, copy_def based on when_def
oheimb
parents: 1461
diff changeset
   126
			   Bound (2*recs_cnt-i) $ Bound (recs_cnt-i);
15574
b1d1b5bfc464 Removed practically all references to Library.foldr.
skalberg
parents: 15570
diff changeset
   127
	val capps = foldr mk_conj (mk_conj(
11531
d038246a62f2 Renamed functions % and %% to avoid clash with syntax for proof terms.
berghofe
parents: 8438
diff changeset
   128
	   Bound(allargs_cnt+1)===mk_cRep_CFun(%%:con,map (bound_arg allvns) vns1),
15574
b1d1b5bfc464 Removed practically all references to Library.foldr.
skalberg
parents: 15570
diff changeset
   129
	   Bound(allargs_cnt+0)===mk_cRep_CFun(%%:con,map (bound_arg allvns) vns2)))
b1d1b5bfc464 Removed practically all references to Library.foldr.
skalberg
parents: 15570
diff changeset
   130
           (mapn rel_app 1 rec_args);
b1d1b5bfc464 Removed practically all references to Library.foldr.
skalberg
parents: 15570
diff changeset
   131
        in foldr mk_ex (Library.foldr mk_conj 
b1d1b5bfc464 Removed practically all references to Library.foldr.
skalberg
parents: 15570
diff changeset
   132
			      (map (defined o Bound) nonlazy_idxs,capps)) allvns end;
1637
b8a8ae2e5de1 Updated: 01-Mar-96 when functional strictified, copy_def based on when_def
oheimb
parents: 1461
diff changeset
   133
      fun one_comp n (_,cons) =mk_all(x_name(n+1),mk_all(x_name(n+1)^"'",mk_imp(
4755
843b5f159c7e added cproj', and therefore extended prj
oheimb
parents: 4122
diff changeset
   134
	 		proj (Bound 2) eqs n $ Bound 1 $ Bound 0,
1637
b8a8ae2e5de1 Updated: 01-Mar-96 when functional strictified, copy_def based on when_def
oheimb
parents: 1461
diff changeset
   135
         		foldr' mk_disj (mk_conj(Bound 1 === UU,Bound 0 === UU)
b8a8ae2e5de1 Updated: 01-Mar-96 when functional strictified, copy_def based on when_def
oheimb
parents: 1461
diff changeset
   136
					::map one_con cons))));
1274
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
   137
    in foldr' mk_conj (mapn one_comp 0 eqs)end ));
16332
25a440fe5f65 add_axioms_infer -- avoids use of stale theory;
wenzelm
parents: 16224
diff changeset
   138
  fun add_one (thy,(dnam,axs,dfs)) = thy
4043
35766855f344 domain package:
oheimb
parents: 4008
diff changeset
   139
	|> Theory.add_path dnam
16332
25a440fe5f65 add_axioms_infer -- avoids use of stale theory;
wenzelm
parents: 16224
diff changeset
   140
	|> add_axioms_infer dfs(*add_defs_i*)
25a440fe5f65 add_axioms_infer -- avoids use of stale theory;
wenzelm
parents: 16224
diff changeset
   141
	|> add_axioms_infer axs
4862
613ce4cc303f adapted to new PureThy.add_axioms_i;
wenzelm
parents: 4755
diff changeset
   142
	|> Theory.parent_path;
15570
8d8c70b41bab Move towards standard functions.
skalberg
parents: 14981
diff changeset
   143
  val thy = Library.foldl add_one (thy', mapn (calc_axioms comp_dname eqs) 0 eqs);
4043
35766855f344 domain package:
oheimb
parents: 4008
diff changeset
   144
in thy |> Theory.add_path comp_dnam  
16332
25a440fe5f65 add_axioms_infer -- avoids use of stale theory;
wenzelm
parents: 16224
diff changeset
   145
       |> add_axioms_infer (bisim_def::(if length eqs>1 then [copy_def] else []))
4862
613ce4cc303f adapted to new PureThy.add_axioms_i;
wenzelm
parents: 4755
diff changeset
   146
       |> Theory.parent_path
4043
35766855f344 domain package:
oheimb
parents: 4008
diff changeset
   147
end;
1274
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
   148
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
   149
end; (* local *)
ea0668a1c0ba added 8bit pragmas
regensbu
parents:
diff changeset
   150
end; (* struct *)