src/HOL/Recdef.thy
author paulson
Tue, 21 Sep 1999 11:11:09 +0200
changeset 7547 a72a551b6d79
parent 7357 d0e16da40ea2
child 7701 2c8c3b7003e5
permissions -rw-r--r--
new proof of drop_prog_correct for new definition of project_act
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
5123
97c1d5c7b701 stepping stones;
wenzelm
parents:
diff changeset
     1
7357
d0e16da40ea2 proper bootstrap of HOL theory and packages;
wenzelm
parents: 6438
diff changeset
     2
theory Recdef = WF_Rel
d0e16da40ea2 proper bootstrap of HOL theory and packages;
wenzelm
parents: 6438
diff changeset
     3
files "Tools/recdef_package.ML" "Tools/induct_method.ML":
6438
e55a1869ed38 'HOL/recdef' theory data;
wenzelm
parents: 5123
diff changeset
     4
e55a1869ed38 'HOL/recdef' theory data;
wenzelm
parents: 5123
diff changeset
     5
setup RecdefPackage.setup
e55a1869ed38 'HOL/recdef' theory data;
wenzelm
parents: 5123
diff changeset
     6
setup InductMethod.setup
e55a1869ed38 'HOL/recdef' theory data;
wenzelm
parents: 5123
diff changeset
     7
e55a1869ed38 'HOL/recdef' theory data;
wenzelm
parents: 5123
diff changeset
     8
end