src/FOL/ex/.if.thy.ML
author nipkow
Mon, 06 Aug 2001 13:43:24 +0200
changeset 11464 ddea204de5bc
parent 0 a5a9c433f639
permissions -rw-r--r--
turned translation for 1::nat into def. introduced 1' and replaced most occurrences of 1 by 1'.

structure If =
struct

local
 val parse_ast_translation = []
 val parse_preproc = None
 val parse_postproc = None
 val parse_translation = []
 val print_translation = []
 val print_preproc = None
 val print_postproc = None
 val print_ast_translation = []
in

(**** begin of user section ****)

(**** end of user section ****)

val thy = extend_theory (FOL.thy)
 "If"
 ([],
  [],
  [],
  [],
  [(["if"], "[o,o,o]=>o")],
  None)
 [("if_def", "if(P,Q,R) == P&Q | ~P&R")]

val ax = get_axiom thy

val if_def = ax "if_def"


end
end